src/HOL/Hilbert_Choice.thy
changeset 58092 4ae52c60603a
parent 58074 87a8cc594bf6
child 58481 62bc7c79212b
--- a/src/HOL/Hilbert_Choice.thy	Thu Aug 28 23:48:46 2014 +0200
+++ b/src/HOL/Hilbert_Choice.thy	Thu Aug 28 23:57:26 2014 +0200
@@ -114,14 +114,14 @@
 subsection {* A skolemization tactic and proof method *}
 
 ML {*
-fun skolem_tac ctxt =
+fun moura_tac ctxt =
   Atomize_Elim.atomize_elim_tac ctxt THEN'
   SELECT_GOAL (Clasimp.auto_tac (ctxt addSIs @{thms choice bchoice}) THEN ALLGOALS (blast_tac ctxt));
 *}
 
-method_setup skolem = {*
- Scan.succeed (SIMPLE_METHOD' o skolem_tac)
-*} "solve skolemization goals"
+method_setup moura = {*
+ Scan.succeed (SIMPLE_METHOD' o moura_tac)
+*} "solve skolemization goals, especially those arising from Z3 proofs"
 
 
 subsection {*Function Inverse*}