# HG changeset patch # User wenzelm # Date 1728395051 -7200 # Node ID 5b201b24d99bec339f336b5c86b751eb4d81b2a9 # Parent 12990a6dddcb01059fc6660e2d97932b79411907 tuned whitespace, to simplify hypersearch; diff -r 12990a6dddcb -r 5b201b24d99b src/Doc/Datatypes/Datatypes.thy --- a/src/Doc/Datatypes/Datatypes.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/Doc/Datatypes/Datatypes.thy Tue Oct 08 15:44:11 2024 +0200 @@ -360,9 +360,7 @@ "[x, xs]" == "x # [xs]" "[x]" == "x # []" - no_notation - Nil (\[]\) and - Cons (infixr \#\ 65) + no_notation Nil (\[]\) and Cons (infixr \#\ 65) hide_type list hide_const Nil Cons case_list hd tl set map list_all2 rec_list size_list list_all diff -r 12990a6dddcb -r 5b201b24d99b src/Doc/Tutorial/ToyList/ToyList.thy --- a/src/Doc/Tutorial/ToyList/ToyList.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/Doc/Tutorial/ToyList/ToyList.thy Tue Oct 08 15:44:11 2024 +0200 @@ -9,7 +9,7 @@ the concrete syntax and name space of theory \<^theory>\Main\ as follows. \ -no_notation Nil ("[]") and Cons (infixr "#" 65) and append (infixr "@" 65) +no_notation Nil ("[]") and Cons (infixr "#" 65) and append (infixr "@" 65) hide_type list hide_const rev diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Analysis/Borel_Space.thy --- a/src/HOL/Analysis/Borel_Space.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Analysis/Borel_Space.thy Tue Oct 08 15:44:11 2024 +0200 @@ -1853,8 +1853,7 @@ shows "f \ borel_measurable M \ g \ borel_measurable M \ Measurable.pred M (\w. f w < g w)" unfolding Measurable.pred_def by (rule borel_measurable_less) -no_notation - eucl_less (infix \ 50) +no_notation eucl_less (infix \ 50) lemma borel_measurable_Max2[measurable (raw)]: fixes f::"_ \ _ \ 'a::{second_countable_topology, dense_linorder, linorder_topology}" diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Analysis/Ordered_Euclidean_Space.thy --- a/src/HOL/Analysis/Ordered_Euclidean_Space.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Analysis/Ordered_Euclidean_Space.thy Tue Oct 08 15:44:11 2024 +0200 @@ -288,8 +288,7 @@ shows "compact {a .. b}" by (metis compact_cbox interval_cbox) -no_notation - eucl_less (infix \ 50) +no_notation eucl_less (infix \ 50) lemma One_nonneg: "0 \ (\Basis::'a::ordered_euclidean_space)" by (auto intro: sum_nonneg) diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Analysis/Topology_Euclidean_Space.thy --- a/src/HOL/Analysis/Topology_Euclidean_Space.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Analysis/Topology_Euclidean_Space.thy Tue Oct 08 15:44:11 2024 +0200 @@ -2484,7 +2484,6 @@ qed qed auto -no_notation - eucl_less (infix \ 50) +no_notation eucl_less (infix \ 50) end diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Examples/Coherent.thy --- a/src/HOL/Examples/Coherent.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Examples/Coherent.thy Tue Oct 08 15:44:11 2024 +0200 @@ -11,9 +11,7 @@ subsection \Equivalence of two versions of Pappus' Axiom\ -no_notation - comp (infixl \o\ 55) and - relcomp (infixr \O\ 75) +no_notation comp (infixl \o\ 55) and relcomp (infixr \O\ 75) lemma p1p2: assumes "col a b c l \ col d e f m" diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Induct/SList.thy --- a/src/HOL/Induct/SList.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Induct/SList.thy Tue Oct 08 15:44:11 2024 +0200 @@ -83,9 +83,7 @@ no_translations "[x, xs]" == "x#[xs]" "[x]" == "x#[]" -no_notation - Nil (\[]\) and - Cons (infixr \#\ 65) +no_notation Nil (\[]\) and Cons (infixr \#\ 65) definition Nil :: "'a list" (\[]\) where diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Library/FSet.thy --- a/src/HOL/Library/FSet.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Library/FSet.thy Tue Oct 08 15:44:11 2024 +0200 @@ -1957,7 +1957,7 @@ end -no_notation Quickcheck_Exhaustive.orelse (infixr \orelse\ 55) +no_notation Quickcheck_Exhaustive.orelse (infixr \orelse\ 55) instantiation fset :: (random) random begin diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Predicate.thy --- a/src/HOL/Predicate.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Predicate.thy Tue Oct 08 15:44:11 2024 +0200 @@ -727,8 +727,7 @@ "pred_of_set (set xs) = foldr sup (List.map Predicate.single xs) bot" by (simp add: pred_of_set_set_fold_sup ac_simps foldr_fold fun_eq_iff) -no_notation - bind (infixl \\\ 70) +no_notation bind (infixl \\\ 70) hide_type (open) pred seq hide_const (open) Pred eval single bind is_empty singleton if_pred not_pred holds diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Probability/ex/Koepf_Duermuth_Countermeasure.thy --- a/src/HOL/Probability/ex/Koepf_Duermuth_Countermeasure.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Probability/ex/Koepf_Duermuth_Countermeasure.thy Tue Oct 08 15:44:11 2024 +0200 @@ -219,7 +219,7 @@ abbreviation joint_probability (\\

'(_ ; _') _\) where "\

(X ; Y) x \ \

(\x. (X x, Y x)) x" -no_notation disj (infixr \|\ 30) +no_notation disj (infixr \|\ 30) abbreviation conditional_probability (\\

'(_ | _') _\) where "\

(X | Y) x \ (\

(X ; Y) x) / \

(Y) (snd`x)" diff -r 12990a6dddcb -r 5b201b24d99b src/HOL/Quotient.thy --- a/src/HOL/Quotient.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/HOL/Quotient.thy Tue Oct 08 15:44:11 2024 +0200 @@ -745,8 +745,7 @@ \Scan.succeed Quotient_Tacs.lifted_attrib\ \lift theorems to quotient types\ -no_notation - rel_conj (infixr \OOO\ 75) +no_notation rel_conj (infixr \OOO\ 75) section \Lifting of BNFs\ diff -r 12990a6dddcb -r 5b201b24d99b src/ZF/ex/Ring.thy --- a/src/ZF/ex/Ring.thy Tue Oct 08 15:02:17 2024 +0200 +++ b/src/ZF/ex/Ring.thy Tue Oct 08 15:44:11 2024 +0200 @@ -6,9 +6,7 @@ theory Ring imports Group begin -no_notation - cadd (infixl \\\ 65) and - cmult (infixl \\\ 70) +no_notation cadd (infixl \\\ 65) and cmult (infixl \\\ 70) (*First, we must simulate a record declaration: record ring = monoid +