This repository has been archived by the owner on Aug 24, 2024. It is now read-only.
-
Notifications
You must be signed in to change notification settings - Fork 16
Commit
This commit does not belong to any branch on this repository, and may belong to a fork outside of the repository.
- Loading branch information
1 parent
de55389
commit 0c4d564
Showing
3 changed files
with
14 additions
and
2 deletions.
There are no files selected for viewing
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1,13 @@ | ||
/-| | ||
Hello World! | ||
-/ | ||
#print "Hello World!" | ||
|
||
/-| | ||
A literate comment! | ||
-/ | ||
|
||
theorem exampleTheorem (p q : Prop) (hp : p) (hq : q) : p ∧ q ∧ p := by | ||
apply And.intro | ||
. exact hp | ||
. sorry |
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1 @@ | ||
[{"contents":[{"typeinfo":null,"semanticType":null,"raw":"/-| \nHello World!\n-/\n","link":null,"docstring":null,"_type":"token"}],"_type":"text"},{"messages":[{"contents":"Hello World!","_type":"message"}],"goals":[],"contents":[{"typeinfo":null,"semanticType":"Keyword","raw":"#print","link":null,"docstring":null,"_type":"token"}],"_type":"sentence"},{"contents":[{"typeinfo":null,"semanticType":null,"raw":" \"Hello World!\"\n\n/-|\nA literate comment!\n-/\n\n","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":"Keyword","raw":"theorem","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" ","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"∀ (p q : Prop), p → q → p ∧ q ∧ p","name":"exampleTheorem","_type":"typeinfo"},"semanticType":null,"raw":"exampleTheorem","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" (","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"Prop","name":"p","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"p","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" ","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"Prop","name":"q","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"q","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" : ","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"Type","name":"Prop","_type":"typeinfo"},"semanticType":null,"raw":"Prop","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":") (","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"p","name":"hp","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"hp","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" : ","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"Prop","name":"p","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"p","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":") (","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"q","name":"hq","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"hq","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" : ","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"Prop","name":"q","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"q","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":") : ","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"Prop","name":"p","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"p","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" ∧ ","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"Prop","name":"q","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"q","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" ∧ ","link":null,"docstring":null,"_type":"token"},{"typeinfo":{"type":"Prop","name":"p","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"p","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" := ","link":null,"docstring":null,"_type":"token"}],"_type":"text"},{"messages":[],"goals":[{"name":"","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"p ∧ q ∧ p","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":"Keyword","raw":"by","link":null,"docstring":null,"_type":"token"},{"typeinfo":null,"semanticType":null,"raw":"\n ","link":null,"docstring":null,"_type":"token"}],"_type":"sentence"},{"messages":[],"goals":[{"name":"left","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"p","_type":"goal"},{"name":"right","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"q ∧ p","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":"Keyword","raw":"apply","link":null,"docstring":"`apply e` tries to match the current goal against the conclusion of `e`'s type.\nIf it succeeds, then the tactic returns as many subgoals as the number of premises that\nhave not been fixed by type inference or type class resolution.\nNon-dependent premises are added before dependent ones.\n\nThe `apply` tactic uses higher-order pattern matching, type class resolution, and first-order unification with dependent types.\n","_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" ","link":null,"docstring":"`apply e` tries to match the current goal against the conclusion of `e`'s type.\nIf it succeeds, then the tactic returns as many subgoals as the number of premises that\nhave not been fixed by type inference or type class resolution.\nNon-dependent premises are added before dependent ones.\n\nThe `apply` tactic uses higher-order pattern matching, type class resolution, and first-order unification with dependent types.\n","_type":"token"},{"typeinfo":{"type":"∀ {a b : Prop}, a → b → a ∧ b","name":"And.intro","_type":"typeinfo"},"semanticType":null,"raw":"And.intro","link":null,"docstring":null,"_type":"token"}],"_type":"sentence"},{"messages":[],"goals":[{"name":"","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"p ∧ q ∧ p","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":null,"raw":"\n ","link":null,"docstring":null,"_type":"token"}],"_type":"sentence"},{"messages":[],"goals":[{"name":"left","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"p","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":null,"raw":".","link":null,"docstring":"`· tac` focuses on the main goal and tries to solve it using `tac`, or else fails. ","_type":"token"}],"_type":"sentence"},{"messages":[],"goals":[{"name":"left","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"p","_type":"goal"},{"name":"right","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"q ∧ p","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":null,"raw":" ","link":null,"docstring":"`· tac` focuses on the main goal and tries to solve it using `tac`, or else fails. ","_type":"token"}],"_type":"sentence"},{"messages":[],"goals":[{"name":"","hypotheses":[],"conclusion":"Goals accomplished! 🐙","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":"Keyword","raw":"exact","link":null,"docstring":"`exact e` closes the main goal if its target type matches that of `e`.\n","_type":"token"},{"typeinfo":null,"semanticType":null,"raw":" ","link":null,"docstring":"`exact e` closes the main goal if its target type matches that of `e`.\n","_type":"token"},{"typeinfo":{"type":"p","name":"hp","_type":"typeinfo"},"semanticType":"Name.Variable","raw":"hp","link":null,"docstring":null,"_type":"token"}],"_type":"sentence"},{"messages":[],"goals":[{"name":"","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"p ∧ q ∧ p","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":null,"raw":"\n ","link":null,"docstring":null,"_type":"token"}],"_type":"sentence"},{"messages":[],"goals":[{"name":"right","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"q ∧ p","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":null,"raw":".","link":null,"docstring":"`· tac` focuses on the main goal and tries to solve it using `tac`, or else fails. ","_type":"token"}],"_type":"sentence"},{"messages":[],"goals":[{"name":"right","hypotheses":[{"type":"Prop","names":["p","q"],"body":"","_type":"hypothesis"},{"type":"p","names":["hp"],"body":"","_type":"hypothesis"},{"type":"q","names":["hq"],"body":"","_type":"hypothesis"}],"conclusion":"q ∧ p","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":null,"raw":" ","link":null,"docstring":"`· tac` focuses on the main goal and tries to solve it using `tac`, or else fails. ","_type":"token"}],"_type":"sentence"},{"messages":[{"contents":"Warning: declaration uses 'sorry'","_type":"message"}],"goals":[{"name":"","hypotheses":[],"conclusion":"Goals accomplished! 🐙","_type":"goal"}],"contents":[{"typeinfo":null,"semanticType":"Keyword","raw":"sorry","link":null,"docstring":"The `sorry` tactic is a shorthand for `exact sorry`. ","_type":"token"}],"_type":"sentence"},{"contents":[],"_type":"text"}] |