src/HOL/Analysis/Simplex_Content.thy
changeset 69173 38beaaebe736
parent 68625 2ec84498f562
child 69517 dc20f278e8f3
--- a/src/HOL/Analysis/Simplex_Content.thy	Sun Oct 21 20:45:01 2018 +0200
+++ b/src/HOL/Analysis/Simplex_Content.thy	Sun Oct 21 23:02:52 2018 +0100
@@ -5,7 +5,7 @@
    The content of an n-dimensional simplex, including the formula for the content of a
    triangle and Heron's formula.
 *)
-section \<open>Volume of a simplex\<close>
+section%important \<open>Volume of a simplex\<close>
 theory Simplex_Content
   imports Change_Of_Vars
 begin
@@ -27,13 +27,13 @@
   using assms sum_nonneg[of A x] unfolding S_def
   by (force simp: sum_delta_notmem algebra_simps)
 
-lemma emeasure_std_simplex_aux:
+lemma%important emeasure_std_simplex_aux:
   fixes t :: real
   assumes "finite (A :: 'a set)" "t \<ge> 0"
   shows   "emeasure (Pi\<^sub>M A (\<lambda>_. lborel)) 
              (S A t \<inter> space (Pi\<^sub>M A (\<lambda>_. lborel))) = t ^ card A / fact (card A)"
   using assms(1,2)
-proof (induction arbitrary: t rule: finite_induct)
+proof%unimportant (induction arbitrary: t rule: finite_induct)
   case (empty t)
   thus ?case by (simp add: PiM_empty S_def)
 next
@@ -111,18 +111,18 @@
   finally show ?thesis by (simp only: std_simplex)
 qed
 
-theorem content_std_simplex:
+theorem%important content_std_simplex:
   "measure lborel (convex hull (insert 0 Basis :: 'a :: euclidean_space set)) =
      1 / fact DIM('a)"
-  by (simp add: measure_def emeasure_std_simplex)
+  by%unimportant (simp add: measure_def emeasure_std_simplex)
 
 (* TODO: move to Change_of_Vars *)
-lemma measure_lebesgue_linear_transformation:
+lemma%important measure_lebesgue_linear_transformation:
   fixes A :: "(real ^ 'n :: {finite, wellorder}) set"
   fixes f :: "_ \<Rightarrow> real ^ 'n :: {finite, wellorder}"
   assumes "bounded A" "A \<in> sets lebesgue" "linear f"
   shows   "measure lebesgue (f ` A) = \<bar>det (matrix f)\<bar> * measure lebesgue A"
-proof -
+proof%unimportant -
   from assms have [intro]: "A \<in> lmeasurable"
     by (intro bounded_set_imp_lmeasurable) auto
   hence [intro]: "f ` A \<in> lmeasurable"
@@ -142,12 +142,12 @@
   finally show ?thesis .
 qed
 
-theorem content_simplex:
+theorem%important content_simplex:
   fixes X :: "(real ^ 'n :: {finite, wellorder}) set" and f :: "'n :: _ \<Rightarrow> real ^ ('n :: _)"
   assumes "finite X" "card X = Suc CARD('n)" and x0: "x0 \<in> X" and bij: "bij_betw f UNIV (X - {x0})"
   defines "M \<equiv> (\<chi> i. \<chi> j. f j $ i - x0 $ i)"
   shows "content (convex hull X) = \<bar>det M\<bar> / fact (CARD('n))"
-proof -
+proof%unimportant -
   define g where "g = (\<lambda>x. M *v x)"
   have [simp]: "M *v axis i 1 = f i - x0" for i :: 'n
     by (simp add: M_def matrix_vector_mult_basis column_def vec_eq_iff)
@@ -183,11 +183,11 @@
     using finite_imp_compact_convex_hull[OF \<open>finite X\<close>] by (auto dest: compact_imp_closed)
 qed
 
-theorem content_triangle:
+theorem%important content_triangle:
   fixes A B C :: "real ^ 2"
   shows "content (convex hull {A, B, C}) =
            \<bar>(C $ 1 - A $ 1) * (B $ 2 - A $ 2) - (B $ 1 - A $ 1) * (C $ 2 - A $ 2)\<bar> / 2"
-proof -
+proof%unimportant -
   define M :: "real ^ 2 ^ 2" where "M \<equiv> (\<chi> i. \<chi> j. (if j = 1 then B else C) $ i - A $ i)"
   define g where "g = (\<lambda>x. M *v x)"
   define std where "std = (convex hull insert 0 Basis :: (real ^ 2) set)"
@@ -227,12 +227,12 @@
     by (auto dest!: compact_imp_closed simp: det_2 M_def)
 qed
 
-theorem heron:
+theorem%important heron:
   fixes A B C :: "real ^ 2"
   defines "a \<equiv> dist B C" and "b \<equiv> dist A C" and "c \<equiv> dist A B"
   defines "s \<equiv> (a + b + c) / 2"
   shows   "content (convex hull {A, B, C}) = sqrt (s * (s - a) * (s - b) * (s - c))"
-proof -
+proof%unimportant -
   have [simp]: "(UNIV :: 2 set) = {1, 2}"
     using exhaust_2 by auto
   have dist_eq: "dist (A :: real ^ 2) B ^ 2 = (A $ 1 - B $ 1) ^ 2 + (A $ 2 - B $ 2) ^ 2"