avoid 'hence' and 'thus' in generated proofs
authorblanchet
Mon, 30 Nov 2015 13:16:12 +0100
changeset 61756 21c2b1f691d1
parent 61755 6af17b2b773d
child 61757 0d399131008f
avoid 'hence' and 'thus' in generated proofs
src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML	Mon Nov 30 13:14:56 2015 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML	Mon Nov 30 13:16:12 2015 +0100
@@ -289,7 +289,7 @@
        else "") ^ "obtain"
 
     fun of_show_have qs = if member (op =) qs Show then "show" else "have"
-    fun of_thus_hence qs = if member (op =) qs Show then "thus" else "hence"
+    fun of_thus_hence qs = if member (op =) qs Show then "then show" else "then have"
 
     fun of_have qs nr =
       if nr > 1 orelse (nr = 1 andalso member (op =) qs Then) then "ultimately " ^ of_show_have qs
@@ -310,8 +310,8 @@
 
     (* Local facts are always passed via "using", which affects "meson" and "metis". This is
        arguably stylistically superior, because it emphasises the structure of the proof. It is also
-       more robust w.r.t. preplay: Preplay is performed before chaining of local facts with "hence"
-       and "thus" is introduced. See also "tac_of_method" in "Sledgehammer_Isar_Preplay". *)
+       more robust w.r.t. preplay: Preplay is performed before chaining of local facts with "then"
+       is introduced. See also "tac_of_method" in "Sledgehammer_Isar_Preplay". *)
     fun of_method ls ss meth =
       let val direct = is_proof_method_direct meth in
         using_facts ls (if direct then [] else ss) ^