# HG changeset patch # User wenzelm # Date 1515359754 -3600 # Node ID 7360fe6bb423acd25202e38745d10aaa47e48db1 # Parent e9bee1ddfe19c1cd5652b25fc35ee4cf72b7f17f prefer formal comments; diff -r e9bee1ddfe19 -r 7360fe6bb423 src/Doc/Isar_Ref/Synopsis.thy --- a/src/Doc/Isar_Ref/Synopsis.thy Sun Jan 07 21:32:21 2018 +0100 +++ b/src/Doc/Isar_Ref/Synopsis.thy Sun Jan 07 22:15:54 2018 +0100 @@ -952,10 +952,10 @@ notepad begin assume r: - "A\<^sub>1 \ A\<^sub>2 \ (* assumptions *) - (\x y. B\<^sub>1 x y \ C\<^sub>1 x y \ R) \ (* case 1 *) - (\x y. B\<^sub>2 x y \ C\<^sub>2 x y \ R) \ (* case 2 *) - R (* main conclusion *)" + "A\<^sub>1 \ A\<^sub>2 \ \ \assumptions\ + (\x y. B\<^sub>1 x y \ C\<^sub>1 x y \ R) \ \ \case 1\ + (\x y. B\<^sub>2 x y \ C\<^sub>2 x y \ R) \ \ \case 2\ + R \ \main conclusion\" have A\<^sub>1 and A\<^sub>2 \ then have R diff -r e9bee1ddfe19 -r 7360fe6bb423 src/HOL/Computational_Algebra/Polynomial.thy --- a/src/HOL/Computational_Algebra/Polynomial.thy Sun Jan 07 21:32:21 2018 +0100 +++ b/src/HOL/Computational_Algebra/Polynomial.thy Sun Jan 07 22:15:54 2018 +0100 @@ -2893,7 +2893,7 @@ where "divide_poly_main lc q r d dr (Suc n) = (let cr = coeff r dr; a = cr div lc; mon = monom a n in - if False \ a * lc = cr then (* False \ is only because of problem in function-package *) + if False \ a * lc = cr then \ \\False \\ is only because of problem in function-package\ divide_poly_main lc (q + mon) diff -r e9bee1ddfe19 -r 7360fe6bb423 src/HOL/Data_Structures/AA_Set.thy --- a/src/HOL/Data_Structures/AA_Set.thy Sun Jan 07 21:32:21 2018 +0100 +++ b/src/HOL/Data_Structures/AA_Set.thy Sun Jan 07 22:15:54 2018 +0100 @@ -29,7 +29,7 @@ fun split :: "'a aa_tree \ 'a aa_tree" where "split (Node lva t1 a (Node lvb t2 b (Node lvc t3 c t4))) = - (if lva = lvb \ lvb = lvc (* lva = lvc suffices *) + (if lva = lvb \ lvb = lvc \ \\lva = lvc\ suffices\ then Node (lva+1) (Node lva t1 a t2) b (Node lva t3 c t4) else Node lva t1 a (Node lvb t2 b (Node lvc t3 c t4)))" | "split t = t" diff -r e9bee1ddfe19 -r 7360fe6bb423 src/HOL/HOLCF/IOA/ABP/Spec.thy --- a/src/HOL/HOLCF/IOA/ABP/Spec.thy Sun Jan 07 21:32:21 2018 +0100 +++ b/src/HOL/HOLCF/IOA/ABP/Spec.thy Sun Jan 07 22:15:54 2018 +0100 @@ -22,7 +22,7 @@ in case fst(snd(tr)) of - Next => t=s | (* Note that there is condition as in Sender *) + Next => t=s | \ \Note that there is condition as in Sender\ S_msg(m) => t = s@[m] | R_msg(m) => s = (m#t) | S_pkt(pkt) => False | diff -r e9bee1ddfe19 -r 7360fe6bb423 src/HOL/Nitpick_Examples/Hotel_Nits.thy --- a/src/HOL/Nitpick_Examples/Hotel_Nits.thy Sun Jan 07 21:32:21 2018 +0100 +++ b/src/HOL/Nitpick_Examples/Hotel_Nits.thy Sun Jan 07 22:15:54 2018 +0100 @@ -44,7 +44,7 @@ "\s \ reach; (k,k') \ cards s g; roomk s r \ {k,k'}\ \ s\isin := (isin s)(r := isin s r \ {g}), roomk := (roomk s)(r := k'), - safe := (safe s)(r := owns s r = Some g \ isin s r = {} (* \ k' = currk s r *) + safe := (safe s)(r := owns s r = Some g \ isin s r = {} \ \\\ k' = currk s r\\ \ safe s r)\ \ reach" | exit_room: "\s \ reach; g \ isin s r\ \ s\isin := (isin s)(r := isin s r - {g})\ \ reach" diff -r e9bee1ddfe19 -r 7360fe6bb423 src/HOL/Quickcheck_Exhaustive.thy --- a/src/HOL/Quickcheck_Exhaustive.thy Sun Jan 07 21:32:21 2018 +0100 +++ b/src/HOL/Quickcheck_Exhaustive.thy Sun Jan 07 22:15:54 2018 +0100 @@ -725,7 +725,7 @@ Some x \ Some x | None \ full_exhaustive_class.full_exhaustive (\(num, t). f (char_of_nat (nat_of_num num), \_ :: unit. Code_Evaluation.App (Code_Evaluation.Const (STR ''String.Char'') TYPEREP(num \ char)) (t ()))) - (min (i - 1) 8) (* generate at most 8 bits *) + (min (i - 1) 8) \ \generate at most 8 bits\ else None)" instance ..