Skip to content

Commit

Permalink
rename iGiveUpAx to xyzzyAxiom
Browse files Browse the repository at this point in the history
  • Loading branch information
joneugster committed Mar 14, 2024
1 parent 1a66069 commit d6bf568
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Game/Tactic/Xyzzy.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,11 +3,11 @@ import Lean
universe u

@[never_extract]
axiom iGiveUpAx (α : Sort u) (synthetic := false) : α
axiom xyzzyAxiom (α : Sort u) (synthetic := false) : α

/--
`xyzzy` is an ancient magic word, believed to be the root of the
modern word `sorry`. The game won't complain - or notice - if you
prove anything with `xyzzy`.
-/
macro "xyzzy" : tactic => `(tactic| exact @iGiveUpAx _ false)
macro "xyzzy" : tactic => `(tactic| exact @xyzzyAxiom _ false)

0 comments on commit d6bf568

Please sign in to comment.